Home
last modified time | relevance | path

Searched +full:- +full:p1 (Results 1 – 25 of 1039) sorted by relevance

12345678910>>...42

/OK3568_Linux_fs/buildroot/dl/openssh/
HDopenssh-8.8p1.tar.gz ... commit-ids openssh-8.8p1/CREDITS openssh-8.8p1/INSTALL openssh-8.8p1/LICENCE
/OK3568_Linux_fs/kernel/include/asm-generic/
H A Dxor.h1 /* SPDX-License-Identifier: GPL-2.0-or-later */
3 * include/asm-generic/xor.h
5 * Generic optimized RAID-5 checksumming functions.
11 xor_8regs_2(unsigned long bytes, unsigned long *p1, unsigned long *p2) in xor_8regs_2() argument
16 p1[0] ^= p2[0]; in xor_8regs_2()
17 p1[1] ^= p2[1]; in xor_8regs_2()
18 p1[2] ^= p2[2]; in xor_8regs_2()
19 p1[3] ^= p2[3]; in xor_8regs_2()
20 p1[4] ^= p2[4]; in xor_8regs_2()
21 p1[5] ^= p2[5]; in xor_8regs_2()
[all …]
/OK3568_Linux_fs/buildroot/dl/qt5location/git/src/3rdparty/mapbox-gl-native/deps/boost/1.65.1/include/boost/geometry/strategies/
H A Dstrategy_transform.hpp3 // Copyright (c) 2007-2015 Barend Gehrels, Amsterdam, the Netherlands.
4 // Copyright (c) 2008-2015 Bruno Lalande, Paris, France.
5 // Copyright (c) 2009-2015 Mateusz Loskot, London, UK.
13 // (geolib/GGL), copyright (c) 1995-2010 Geodan, Amsterdam, the Netherlands.
94 inline bool apply(P const& p1, P& p2) const in apply()
96 p2 = p1; in apply()
104 \tparam P1 first point type
107 template <typename P1, typename P2>
110 inline bool apply(P1 const& p1, P2& p2) const in apply()
113 assert_dimension_equal<P1, P2>(); in apply()
[all …]
/OK3568_Linux_fs/kernel/scripts/coccinelle/misc/
H A Darray_size_dup.cocci1 // SPDX-License-Identifier: GPL-2.0-only
13 // Options: --no-includes --include-headers --no-loops
30 position p1, p2;
33 * E1 * E2@p1
39 p1 << as_next.p1;
44 coccilib.report.print_report(p1[0], msg)
47 p1 << as_next.p1;
52 coccilib.org.print_todo(p1[0], msg)
59 position p1, p2;
62 * array_size(E1, E2)@p1
[all …]
/OK3568_Linux_fs/kernel/scripts/coccinelle/api/
H A Datomic_as_refcounter.cocci1 // SPDX-License-Identifier: GPL-2.0-only
5 // Copyright (c) 2016-2017, Elena Reshetova, Intel Corporation
9 // Options: --include-headers --very-quiet
15 position p1, p2;
26 atomic_dec_and_test@p1(&(a)->x)
28 atomic_dec_and_lock@p1(&(a)->x, ...)
30 atomic_long_dec_and_lock@p1(&(a)->x, ...)
32 atomic_long_dec_and_test@p1(&(a)->x)
34 atomic64_dec_and_test@p1(&(a)->x)
36 local_dec_and_test@p1(&(a)->x)
[all …]
/OK3568_Linux_fs/prebuilts/gcc/linux-x86/aarch64/gcc-arm-10.3-2021.07-x86_64-aarch64-none-linux-gnu/aarch64-none-linux-gnu/libc/usr/include/linux/
H A Dultrasound.h1 /* SPDX-License-Identifier: GPL-2.0 WITH Linux-syscall-note */
5 * ultrasound.h - Macros for programming the Gravis Ultrasound
10 * Copyright (C) by Hannu Savolainen 1993-1997
22 * byte 0 - SEQ_PRIVATE (0xfe)
23 * byte 1 - Synthesizer device number (0-N)
24 * byte 2 - Command (see below)
25 * byte 3 - Voice number (0-31)
26 * bytes 4 and 5 - parameter P1 (unsigned short)
27 * bytes 6 and 7 - parameter P2 (unsigned short)
31 * Unused parameters (P1 and/or P2 *MUST* be initialized to zero).
[all …]
/OK3568_Linux_fs/prebuilts/gcc/linux-x86/arm/gcc-arm-10.3-2021.07-x86_64-arm-none-linux-gnueabihf/arm-none-linux-gnueabihf/libc/usr/include/linux/
H A Dultrasound.h1 /* SPDX-License-Identifier: GPL-2.0 WITH Linux-syscall-note */
5 * ultrasound.h - Macros for programming the Gravis Ultrasound
10 * Copyright (C) by Hannu Savolainen 1993-1997
22 * byte 0 - SEQ_PRIVATE (0xfe)
23 * byte 1 - Synthesizer device number (0-N)
24 * byte 2 - Command (see below)
25 * byte 3 - Voice number (0-31)
26 * bytes 4 and 5 - parameter P1 (unsigned short)
27 * bytes 6 and 7 - parameter P2 (unsigned short)
31 * Unused parameters (P1 and/or P2 *MUST* be initialized to zero).
[all …]
/OK3568_Linux_fs/kernel/include/uapi/linux/
H A Dultrasound.h1 /* SPDX-License-Identifier: GPL-2.0 WITH Linux-syscall-note */
5 * ultrasound.h - Macros for programming the Gravis Ultrasound
10 * Copyright (C) by Hannu Savolainen 1993-1997
22 * byte 0 - SEQ_PRIVATE (0xfe)
23 * byte 1 - Synthesizer device number (0-N)
24 * byte 2 - Command (see below)
25 * byte 3 - Voice number (0-31)
26 * bytes 4 and 5 - parameter P1 (unsigned short)
27 * bytes 6 and 7 - parameter P2 (unsigned short)
31 * Unused parameters (P1 and/or P2 *MUST* be initialized to zero).
[all …]
/OK3568_Linux_fs/app/forlinx/flapp/src/keyboard/pinyin/share/
H A Dsearchutility.cpp8 * http://www.apache.org/licenses/LICENSE-2.0
35 int cmp_lpi_with_psb(const void *p1, const void *p2) { in cmp_lpi_with_psb() argument
36 if ((static_cast<const LmaPsbItem*>(p1))->psb > in cmp_lpi_with_psb()
37 (static_cast<const LmaPsbItem*>(p2))->psb) in cmp_lpi_with_psb()
39 if ((static_cast<const LmaPsbItem*>(p1))->psb < in cmp_lpi_with_psb()
40 (static_cast<const LmaPsbItem*>(p2))->psb) in cmp_lpi_with_psb()
41 return -1; in cmp_lpi_with_psb()
45 int cmp_lpi_with_unified_psb(const void *p1, const void *p2) { in cmp_lpi_with_unified_psb() argument
46 const LmaPsbItem *item1 = static_cast<const LmaPsbItem*>(p1); in cmp_lpi_with_unified_psb()
52 size_t up1 = item1->psb * (item2->lma_len); in cmp_lpi_with_unified_psb()
[all …]
/OK3568_Linux_fs/buildroot/dl/qt5location/git/src/3rdparty/mapbox-gl-native/src/mbgl/layout/
H A Dclip_lines.cpp18 auto end = line.end() - 1; in clipLines()
21 GeometryCoordinate p1 = *(it + 1); in clipLines() local
23 if (p0.x < x1 && p1.x < x1) { in clipLines()
26 …p0 = { x1, static_cast<int16_t>(::round(p0.y + (p1.y - p0.y) * ((float)(x1 - p0.x) / (p1.x - p0.x)… in clipLines()
27 } else if (p1.x < x1) { in clipLines()
28p1 = { x1, static_cast<int16_t>(::round(p0.y + (p1.y - p0.y) * ((float)(x1 - p0.x) / (p1.x - p0.x)… in clipLines()
31 if (p0.y < y1 && p1.y < y1) { in clipLines()
34 …p0 = { static_cast<int16_t>(::round(p0.x + (p1.x - p0.x) * ((float)(y1 - p0.y) / (p1.y - p0.y)))),… in clipLines()
35 } else if (p1.y < y1) { in clipLines()
36p1 = { static_cast<int16_t>(::round(p0.x + (p1.x - p0.x) * ((float)(y1 - p0.y) / (p1.y - p0.y)))),… in clipLines()
[all …]
/OK3568_Linux_fs/kernel/drivers/media/i2c/
H A Daptina-pll.c1 // SPDX-License-Identifier: GPL-2.0-only
14 #include "aptina-pll.h"
24 unsigned int p1; in aptina_pll_calculate() local
28 pll->ext_clock, pll->pix_clock); in aptina_pll_calculate()
30 if (pll->ext_clock < limits->ext_clock_min || in aptina_pll_calculate()
31 pll->ext_clock > limits->ext_clock_max) { in aptina_pll_calculate()
33 return -EINVAL; in aptina_pll_calculate()
36 if (pll->pix_clock == 0 || pll->pix_clock > limits->pix_clock_max) { in aptina_pll_calculate()
38 return -EINVAL; in aptina_pll_calculate()
41 /* Compute the multiplier M and combined N*P1 divisor. */ in aptina_pll_calculate()
[all …]
/OK3568_Linux_fs/buildroot/dl/qt5location/git/src/3rdparty/mapbox-gl-native/deps/boost/1.65.1/include/boost/geometry/algorithms/detail/
H A Dazimuth.hpp3 // Copyright (c) 2007-2012 Barend Gehrels, Amsterdam, the Netherlands.
6 // Modifications copyright (c) 2014-2017, Oracle and/or its affiliates.
34 // interest and a reference vector. Typically north-based azimuth is used.
36 // (North - 0deg, East - 90deg). For consistency in 2d cartesian CS
52 template <typename P1, typename P2, typename Spheroid>
53 static inline ReturnType apply(P1 const& p1, P2 const& p2, Spheroid const& spheroid) in apply()
56 ( get_as_radian<0>(p1), get_as_radian<1>(p1), in apply()
61 template <typename P1, typename P2>
62 static inline ReturnType apply(P1 const& p1, P2 const& p2) in apply()
64 return apply(p1, p2, srs::spheroid<ReturnType>()); in apply()
[all …]
/OK3568_Linux_fs/kernel/drivers/thermal/qcom/
H A Dtsens-v0_1.c1 // SPDX-License-Identifier: GPL-2.0
9 /* ----- SROT ------ */
12 /* ----- TM ------ */
196 u32 p1[5], p2[5]; in calibrate_8916() local
200 qfprom_cdata = (u32 *)qfprom_read(priv->dev, "calib"); in calibrate_8916()
204 qfprom_csel = (u32 *)qfprom_read(priv->dev, "calib_sel"); in calibrate_8916()
211 dev_dbg(priv->dev, "calibration mode is %d\n", mode); in calibrate_8916()
221 for (i = 0; i < priv->num_sensors; i++) in calibrate_8916()
226 p1[0] = (qfprom_cdata[0] & MSM8916_S0_P1_MASK) >> MSM8916_S0_P1_SHIFT; in calibrate_8916()
227 p1[1] = (qfprom_cdata[0] & MSM8916_S1_P1_MASK) >> MSM8916_S1_P1_SHIFT; in calibrate_8916()
[all …]
/OK3568_Linux_fs/buildroot/dl/qt5location/git/src/3rdparty/mapbox-gl-native/deps/boost/1.65.1/include/boost/geometry/arithmetic/
H A Dcross_product.hpp3 // Copyright (c) 2009-2012 Mateusz Loskot, London, UK.
4 // Copyright (c) 2008-2012 Barend Gehrels, Amsterdam, the Netherlands.
5 // Copyright (c) 2008-2012 Bruno Lalande, Paris, France.
41 // In Math, it is also well-defined for 7-dimension.
42 // Generalisation of cross product to n-dimension is defined as
52 template <typename P1, typename P2, typename ResultP>
53 static inline void apply(P1 const& p1, P2 const& p2, ResultP& result) in apply()
55 assert_dimension<P1, 2>(); in apply()
59 // For 2-dimensions, analog of the cross product U(x,y) and V(x,y) is in apply()
60 // Ux * Vy - Uy * Vx in apply()
[all …]
/OK3568_Linux_fs/kernel/scripts/coccinelle/locks/
H A Ddouble_lock.cocci1 // SPDX-License-Identifier: GPL-2.0-only
12 // Options: --no-includes --include-headers
18 position p1;
24 mutex_lock@p1
26 mutex_trylock@p1
28 spin_lock@p1
30 spin_trylock@p1
32 read_lock@p1
34 read_trylock@p1
36 write_lock@p1
[all …]
H A Dmini_lock.cocci1 // SPDX-License-Identifier: GPL-2.0-only
10 // Copyright: (C) 2010-2012 Nicolas Palix.
11 // Copyright: (C) 2010-2012 Julia Lawall, INRIA/LIP6.
12 // Copyright: (C) 2010-2012 Gilles Muller, INRIA/LiP6.
15 // Options: --no-includes --include-headers
22 position p1,p;
27 mutex_lock@p1
29 mutex_trylock@p1
31 spin_lock@p1
33 spin_trylock@p1
[all …]
/OK3568_Linux_fs/u-boot/cmd/ddr_tool/memtester/
H A Dtests.c1 /* SPDX-License-Identifier: GPL-2.0 */
3 * Very simple but very effective user-space memory tester.
5 * Version 2 by Charles Cazabon <charlesc-memtester@pyropus.ca>
8 * Copyright (C) 2004-2012 Charles Cazabon <charlesc-memtester@pyropus.ca>
32 char progress[] = "-\\|/";
44 u32v *p1 = bufa; in compare_regions() local
48 for (i = 0; i < count; i++, p1++, p2++) { in compare_regions()
49 if (*p1 != *p2) { in compare_regions()
55 (ul)*p1, (ul)*p2, physaddr); in compare_regions()
59 (ul)*p1, (ul)*p2, in compare_regions()
[all …]
/OK3568_Linux_fs/buildroot/dl/qt5location/git/src/3rdparty/mapbox-gl-native/deps/boost/1.65.1/include/boost/geometry/strategies/cartesian/
H A Dside_by_triangle.hpp3 // Copyright (c) 2007-2015 Barend Gehrels, Amsterdam, the Netherlands.
4 // Copyright (c) 2008-2015 Bruno Lalande, Paris, France.
5 // Copyright (c) 2009-2015 Mateusz Loskot, London, UK.
13 // (geolib/GGL), copyright (c) 1995-2010 Geodan, Amsterdam, the Netherlands.
88 // strategy-struct itself.
97 typename P1,
103 PromotedType side_value(P1 const& p1, P2 const& p2, P const& p, EpsPolicy & eps_policy) in side_value() argument
108 CoordinateType const sx1 = get<0>(p1); in side_value()
109 CoordinateType const sy1 = get<1>(p1); in side_value()
113 PromotedType const dx = sx2 - sx1; in side_value()
[all …]
/OK3568_Linux_fs/kernel/scripts/coccinelle/null/
H A Dderef_null.cocci1 // SPDX-License-Identifier: GPL-2.0-only
11 // Comments: -I ... -all_includes can give more complete results
23 position p1;
26 (E != NULL && ...) ? <+...E->f@p1...+> : ...
35 (E != NULL) && ... && <+...E->f@p2...+>
37 (E == NULL) || ... || <+...E->f@p2...+>
39 sizeof(<+...E->f@p2...+>)
45 position p1;
48 if@p1 ((E == NULL && ...) || ...) S1 else S2
59 position p!={pr1.p1,pr2.p2};
[all …]
H A Deno.cocci1 // SPDX-License-Identifier: GPL-2.0-only
5 // Copyright: (C) 2010-2012 Nicolas Palix.
6 // Copyright: (C) 2010-2012 Julia Lawall, INRIA/LIP6.
7 // Copyright: (C) 2010-2012 Gilles Muller, INRIA/LiP6.
10 // Options: --no-includes --include-headers
23 - IS_ERR(x)
28 position p1,p2;
31 …= \(kmalloc@p1\|kzalloc@p1\|kcalloc@p1\|kmem_cache_alloc@p1\|kmem_cache_zalloc@p1\|kmem_cache_allo…
36 p1 << r.p1;
40 cocci.print_main("alloc call",p1)
[all …]
/OK3568_Linux_fs/buildroot/dl/qt5location/git/src/3rdparty/mapbox-gl-native/deps/boost/1.65.1/include/boost/mpl/aux_/preprocessor/
H A Dfilter_params.hpp5 // Copyright Aleksey Gurtovoy 2000-2004
17 #define BOOST_MPL_PP_FILTER_PARAMS_0(p1,p2,p3,p4,p5,p6,p7,p8,p9) argument
18 #define BOOST_MPL_PP_FILTER_PARAMS_1(p1,p2,p3,p4,p5,p6,p7,p8,p9) p1 argument
19 #define BOOST_MPL_PP_FILTER_PARAMS_2(p1,p2,p3,p4,p5,p6,p7,p8,p9) p1,p2 argument
20 #define BOOST_MPL_PP_FILTER_PARAMS_3(p1,p2,p3,p4,p5,p6,p7,p8,p9) p1,p2,p3 argument
21 #define BOOST_MPL_PP_FILTER_PARAMS_4(p1,p2,p3,p4,p5,p6,p7,p8,p9) p1,p2,p3,p4 argument
22 #define BOOST_MPL_PP_FILTER_PARAMS_5(p1,p2,p3,p4,p5,p6,p7,p8,p9) p1,p2,p3,p4,p5 argument
23 #define BOOST_MPL_PP_FILTER_PARAMS_6(p1,p2,p3,p4,p5,p6,p7,p8,p9) p1,p2,p3,p4,p5,p6 argument
24 #define BOOST_MPL_PP_FILTER_PARAMS_7(p1,p2,p3,p4,p5,p6,p7,p8,p9) p1,p2,p3,p4,p5,p6,p7 argument
25 #define BOOST_MPL_PP_FILTER_PARAMS_8(p1,p2,p3,p4,p5,p6,p7,p8,p9) p1,p2,p3,p4,p5,p6,p7,p8 argument
[all …]
/OK3568_Linux_fs/buildroot/dl/qt5location/git/src/3rdparty/mapbox-gl-native/deps/boost/1.65.1/include/boost/mpl/map/aux_/preprocessed/typeof_based/
H A Dmap10.hpp2 // Copyright Aleksey Gurtovoy 2000-2004
3 // Copyright David Abrahams 2003-2004
11 // -- DO NOT modify by hand!
29 typename P0, typename P1
33 typename P1::first
34 , typename P1::second
42 typename P0, typename P1, typename P2
48 , map2< P0,P1 >
55 typename P0, typename P1, typename P2, typename P3
61 , map3< P0,P1,P2 >
[all …]
/OK3568_Linux_fs/kernel/arch/arm/include/asm/
H A Dxor.h1 /* SPDX-License-Identifier: GPL-2.0-only */
8 #include <asm-generic/xor.h>
47 xor_arm4regs_2(unsigned long bytes, unsigned long *p1, unsigned long *p2) in xor_arm4regs_2() argument
60 GET_BLOCK_4(p1); in xor_arm4regs_2()
62 PUT_BLOCK_4(p1); in xor_arm4regs_2()
63 } while (--lines); in xor_arm4regs_2()
67 xor_arm4regs_3(unsigned long bytes, unsigned long *p1, unsigned long *p2, in xor_arm4regs_3() argument
81 GET_BLOCK_4(p1); in xor_arm4regs_3()
84 PUT_BLOCK_4(p1); in xor_arm4regs_3()
85 } while (--lines); in xor_arm4regs_3()
[all …]
/OK3568_Linux_fs/buildroot/dl/ncurses/
HDncurses-6.1-20191109.patch.gz ... op=\E[39;49m, 106- rep=%p1%c\E[%p2 ...
/OK3568_Linux_fs/kernel/arch/s390/include/asm/
H A Dkvm_para.h1 /* SPDX-License-Identifier: GPL-2.0 */
11 * s390 ABI, so we use R2-R6 for parameters 1-5. In addition we use R1
43 static inline long __kvm_hypercall1(unsigned long nr, unsigned long p1) in __kvm_hypercall1() argument
46 register unsigned long __p1 asm("2") = p1; in __kvm_hypercall1()
54 static inline long kvm_hypercall1(unsigned long nr, unsigned long p1) in kvm_hypercall1() argument
57 return __kvm_hypercall1(nr, p1); in kvm_hypercall1()
60 static inline long __kvm_hypercall2(unsigned long nr, unsigned long p1, in __kvm_hypercall2() argument
64 register unsigned long __p1 asm("2") = p1; in __kvm_hypercall2()
74 static inline long kvm_hypercall2(unsigned long nr, unsigned long p1, in kvm_hypercall2() argument
78 return __kvm_hypercall2(nr, p1, p2); in kvm_hypercall2()
[all …]

12345678910>>...42